blob: edecee79e7e5c670ca7e66f5dc5117553a0963fe (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
|
(* Test of inference of elimination predicate for "if" *)
(* submitted by Robert R Schneck *)
Axiom bad : false = true.
Definition try1 : False :=
<[b:bool][_:false=b](if b then False else True)>
Cases bad of refl_equal => I end.
Definition try2 : False :=
<[b:bool][_:false=b]((if b then False else True)::Prop)>
Cases bad of refl_equal => I end.
Definition try3 : False :=
<[b:bool][_:false=b](([b':bool] if b' then False else True) b)>
Cases bad of refl_equal => I end.
|