File: simpl_done.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 (28 lines) | stat: -rw-r--r-- 547 bytes parent folder | download | duplicates (5)
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
Require Import ssreflect.

Inductive lit : Set :=
| LitP : lit
| LitL : lit
.

Inductive val : Set :=
| Val : lit -> val.

Definition tyref :=
fun (vl : list val) =>
match vl with
| cons (Val LitL) (cons (Val LitP) _)  => False
| _ => False
end.

(** Check that simplification and resolution are performed in the right order
    by "//=" when several goals are under focus. *)
Goal exists vl1 : list val,
  cons (Val LitL) (cons (Val LitL) nil) = vl1 /\
  (tyref vl1)
.
Proof.
eexists (cons _ (cons _ _)).
split =>//=.
Fail progress simpl.
Abort.