File: bug_18503.v

package info (click to toggle)
coq 8.20.1%2Bdfsg-1
  • links: PTS, VCS
  • area: main
  • in suites: sid, trixie
  • size: 44,116 kB
  • sloc: ml: 234,160; sh: 4,301; python: 3,270; ansic: 2,644; makefile: 882; lisp: 172; javascript: 63; xml: 24; sed: 2
file content (41 lines) | stat: -rw-r--r-- 659 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
Require Import PrimInt63.
Open Scope int63_scope.

Module Type T.
  Primitive bar := #int63_sub.

  Axiom bar_land : bar = land.
End T.

Module F(X:T).
  Definition foo : X.bar 1 1 = 0 := eq_refl.
End F.

Module M.
  Definition bar := land.
  Definition bar_land : bar = land := eq_refl.
End M.

Fail Module N : T := M.

(*
Module A := F N.

Lemma bad : False.
Proof.
  pose (f := fun x => eqb x 1).
  assert (H:f 1 = f 0).
  { f_equal. change 1 with (land 1 1).
    rewrite <-N.bar_land.
    exact A.foo. }
  change (true = false) in H.
  inversion H.
Qed.

Print Assumptions bad.
(* Axioms:
land : int -> int -> int
int : Set
eqb : int -> int -> bool
*)
*)