Nominal/Term5.thy
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Sat, 20 Mar 2010 10:12:09 +0100
changeset 1562 41294e4fc870
parent 1489 b9caceeec805
child 1575 2c37f5a8c747
permissions -rw-r--r--
Size experiments.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     1
theory Term5
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     2
imports "Nominal2_Atoms" "Nominal2_Eqvt" "Nominal2_Supp" "Abs" "Perm" "Fv" "Rsp" "../Attic/Prove"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     3
begin
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     4
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     5
atom_decl name
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     6
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     7
datatype rtrm5 =
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     8
  rVr5 "name"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
     9
| rAp5 "rtrm5" "rtrm5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    10
| rLt5 "rlts" "rtrm5" --"bind (bv5 lts) in (rtrm5)"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    11
and rlts =
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    12
  rLnil
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    13
| rLcons "name" "rtrm5" "rlts"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    14
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    15
primrec
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    16
  rbv5
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    17
where
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    18
  "rbv5 rLnil = {}"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    19
| "rbv5 (rLcons n t ltl) = {atom n} \<union> (rbv5 ltl)"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    20
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    21
1277
6eacf60ce41d Permutation and FV_Alpha interface change.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1270
diff changeset
    22
setup {* snd o define_raw_perms (Datatype.the_info @{theory} "Term5.rtrm5") 2 *}
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    23
print_theorems
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    24
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
    25
local_setup {* snd o define_fv_alpha (Datatype.the_info @{theory} "Term5.rtrm5")
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
    26
  [[[], [], [(SOME (@{term rbv5}, true), 0, 1)]], [[], []]] [(@{term rbv5}, 1, [[], [0, 2]])] *}
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    27
print_theorems
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    28
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    29
notation
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    30
  alpha_rtrm5 ("_ \<approx>5 _" [100, 100] 100) and
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    31
  alpha_rlts ("_ \<approx>l _" [100, 100] 100)
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
    32
thm alpha_rtrm5_alpha_rlts_alpha_rbv5.intros
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    33
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
    34
local_setup {* (fn ctxt => snd (Local_Theory.note ((@{binding alpha5_inj}, []), (build_alpha_inj @{thms alpha_rtrm5_alpha_rlts_alpha_rbv5.intros} @{thms rtrm5.distinct rtrm5.inject rlts.distinct rlts.inject} @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} ctxt)) ctxt)) *}
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    35
thm alpha5_inj
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    36
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    37
lemma rbv5_eqvt[eqvt]:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    38
  "pi \<bullet> (rbv5 x) = rbv5 (pi \<bullet> x)"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    39
  apply (induct x)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    40
  apply (simp_all add: eqvts atom_eqvt)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    41
  done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    42
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    43
lemma fv_rtrm5_rlts_eqvt[eqvt]:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    44
  "pi \<bullet> (fv_rtrm5 x) = fv_rtrm5 (pi \<bullet> x)"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    45
  "pi \<bullet> (fv_rlts l) = fv_rlts (pi \<bullet> l)"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    46
  apply (induct x and l)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    47
  apply (simp_all add: eqvts atom_eqvt)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    48
  done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    49
1455
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    50
(*lemma alpha5_eqvt:
1419
3cf30bb8c6f6 The alpha5_eqvt tactic works if I manage to build the goal.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1405
diff changeset
    51
  "(xa \<approx>5 y \<longrightarrow> (p \<bullet> xa) \<approx>5 (p \<bullet> y)) \<and>
3cf30bb8c6f6 The alpha5_eqvt tactic works if I manage to build the goal.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1405
diff changeset
    52
  (xb \<approx>l ya \<longrightarrow> (p \<bullet> xb) \<approx>l (p \<bullet> ya)) \<and>
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    53
  (alpha_rbv5 b c \<longrightarrow> alpha_rbv5 (p \<bullet> b) (p \<bullet> c))"
1419
3cf30bb8c6f6 The alpha5_eqvt tactic works if I manage to build the goal.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1405
diff changeset
    54
apply (tactic {* alpha_eqvt_tac @{thm alpha_rtrm5_alpha_rlts_alpha_rbv5.induct} @{thms alpha5_inj permute_rtrm5_permute_rlts.simps} @{context} 1 *})
1455
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    55
done*)
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    56
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    57
local_setup {*
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    58
(fn ctxt => snd (Local_Theory.note ((@{binding alpha5_eqvt}, []),
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    59
build_alpha_eqvts [@{term alpha_rtrm5}, @{term alpha_rlts}, @{term alpha_rbv5}] (fn _ => alpha_eqvt_tac  @{thm alpha_rtrm5_alpha_rlts_alpha_rbv5.induct} @{thms alpha5_inj permute_rtrm5_permute_rlts.simps} ctxt 1) ctxt) ctxt)) *}
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    60
print_theorems
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
    61
1421
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    62
lemma alpha5_reflp:
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
    63
"y \<approx>5 y \<and> (x \<approx>l x \<and> alpha_rbv5 x x)"
1421
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    64
apply (rule rtrm5_rlts.induct)
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    65
apply (simp_all add: alpha5_inj)
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    66
apply (rule_tac x="0::perm" in exI)
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    67
apply (simp add: eqvts alpha_gen fresh_star_def fresh_zero_perm)
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    68
done
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    69
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    70
lemma alpha5_symp:
1453
49bdb8d475df The proof in 'Test' gets simpler.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1421
diff changeset
    71
"(a \<approx>5 b \<longrightarrow> b \<approx>5 a) \<and>
1421
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    72
(x \<approx>l y \<longrightarrow> y \<approx>l x) \<and>
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
    73
(alpha_rbv5 x y \<longrightarrow> alpha_rbv5 y x)"
1489
b9caceeec805 compose_sym2 works also for term5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1474
diff changeset
    74
apply (tactic {* symp_tac @{thm alpha_rtrm5_alpha_rlts_alpha_rbv5.induct} @{thms alpha5_inj} @{thms alpha5_eqvt} @{context} 1 *})
b9caceeec805 compose_sym2 works also for term5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1474
diff changeset
    75
(*
1421
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    76
apply (rule alpha_rtrm5_alpha_rlts_alpha_rbv5.induct)
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
    77
apply (simp_all add: alpha5_inj)
1455
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    78
apply (erule exE)
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    79
apply (rule_tac x="- pi" in exI)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    80
apply (simp add: alpha_gen)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    81
  apply(simp add: fresh_star_def fresh_minus_perm)
1455
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    82
apply clarify
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
    83
apply (rule conjI)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    84
apply (rotate_tac 3)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    85
apply (frule_tac p="- pi" in alpha5_eqvt(2))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    86
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    87
apply (rule conjI)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    88
apply (rotate_tac 5)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    89
apply (frule_tac p="- pi" in alpha5_eqvt(1))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    90
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    91
apply (rotate_tac 6)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    92
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
    93
apply (drule_tac p1="- pi" in permute_eq_iff[symmetric,THEN iffD1])
1489
b9caceeec805 compose_sym2 works also for term5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1474
diff changeset
    94
apply (simp)*)
1455
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    95
done
0fae5608cd1e alpha5_symp proved.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1454
diff changeset
    96
1456
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
    97
lemma alpha5_transp:
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
    98
"(a \<approx>5 b \<longrightarrow> (\<forall>c. b \<approx>5 c \<longrightarrow> a \<approx>5 c)) \<and>
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
    99
(x \<approx>l y \<longrightarrow> (\<forall>z. y \<approx>l z \<longrightarrow> x \<approx>l z)) \<and>
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   100
(alpha_rbv5 k l \<longrightarrow> (\<forall>m. alpha_rbv5 l m \<longrightarrow> alpha_rbv5 k m))"
1456
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   101
(*apply (tactic {* transp_tac @{context} @{thm alpha_rtrm5_alpha_rlts_alpha_rbv5.induct} @{thms alpha5_inj} @{thms rtrm5.distinct rtrm5.inject rlts.distinct rlts.inject} [] @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{thms alpha5_eqvt} 1 *})*)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   102
apply (rule alpha_rtrm5_alpha_rlts_alpha_rbv5.induct)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   103
apply (rule_tac [!] allI)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   104
apply (tactic {* (imp_elim_tac @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{context}) 1 *})
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   105
apply (simp_all add: alpha5_inj)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   106
apply (tactic {* (imp_elim_tac @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{context}) 1 *})
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   107
apply (simp_all add: alpha5_inj)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   108
apply (tactic {* (imp_elim_tac @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{context}) 1 *})
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   109
apply (simp_all add: alpha5_inj)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   110
defer
1456
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   111
apply (tactic {* (imp_elim_tac @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{context}) 1 *})
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   112
apply (simp_all add: alpha5_inj)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   113
apply (tactic {* (imp_elim_tac @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases} @{context}) 1 *})
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   114
apply (simp_all add: alpha5_inj)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   115
apply (tactic {* eetac @{thm exi_sum} @{context} 1 *})
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   116
apply (simp add: alpha_gen)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   117
apply clarify
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   118
apply(simp add: fresh_star_plus)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   119
apply (rule conjI)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   120
apply (erule_tac x="- pi \<bullet> rltsaa" in allE)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   121
apply (rotate_tac 5)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   122
apply (drule_tac p="- pi" in alpha5_eqvt(2))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   123
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   124
apply (drule_tac p="pi" in alpha5_eqvt(2))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   125
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   126
apply (erule_tac x="- pi \<bullet> rtrm5aa" in allE)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   127
apply (rotate_tac 7)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   128
apply (drule_tac p="- pi" in alpha5_eqvt(1))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   129
apply simp
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   130
apply (rotate_tac 3)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   131
apply (drule_tac p="pi" in alpha5_eqvt(1))
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   132
apply simp
1456
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   133
done
1421
95324fb345e5 looking at trm5_equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1419
diff changeset
   134
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   135
lemma alpha5_equivp:
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   136
  "equivp alpha_rtrm5"
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   137
  "equivp alpha_rlts"
1456
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   138
  unfolding equivp_reflp_symp_transp reflp_def symp_def transp_def
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   139
  apply (simp_all only: alpha5_reflp)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   140
  apply (meson alpha5_symp alpha5_transp)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   141
  apply (meson alpha5_symp alpha5_transp)
686c58ea7a24 alpha5_transp and equivp
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1455
diff changeset
   142
  done
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   143
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   144
quotient_type
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   145
  trm5 = rtrm5 / alpha_rtrm5
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   146
and
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   147
  lts = rlts / alpha_rlts
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   148
  by (auto intro: alpha5_equivp)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   149
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   150
local_setup {*
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   151
(fn ctxt => ctxt
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   152
 |> snd o (Quotient_Def.quotient_lift_const ("Vr5", @{term rVr5}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   153
 |> snd o (Quotient_Def.quotient_lift_const ("Ap5", @{term rAp5}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   154
 |> snd o (Quotient_Def.quotient_lift_const ("Lt5", @{term rLt5}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   155
 |> snd o (Quotient_Def.quotient_lift_const ("Lnil", @{term rLnil}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   156
 |> snd o (Quotient_Def.quotient_lift_const ("Lcons", @{term rLcons}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   157
 |> snd o (Quotient_Def.quotient_lift_const ("fv_trm5", @{term fv_rtrm5}))
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   158
 |> snd o (Quotient_Def.quotient_lift_const ("fv_lts", @{term fv_rlts}))
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   159
 |> snd o (Quotient_Def.quotient_lift_const ("bv5", @{term rbv5}))
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   160
 |> snd o (Quotient_Def.quotient_lift_const ("alpha_bv5", @{term alpha_rbv5})))
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   161
*}
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   162
print_theorems
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   163
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   164
lemma alpha5_rfv:
1405
3e128904baba More tries about the proofs in trm5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1402
diff changeset
   165
  "(t \<approx>5 s \<Longrightarrow> fv_rtrm5 t = fv_rtrm5 s)"
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   166
  "(l \<approx>l m \<Longrightarrow> fv_rlts l = fv_rlts m)"
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   167
  "(alpha_rbv5 b c \<Longrightarrow> True)"
1405
3e128904baba More tries about the proofs in trm5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1402
diff changeset
   168
  apply(induct rule: alpha_rtrm5_alpha_rlts_alpha_rbv5.inducts)
1454
7c8cd6eae8e2 FV_bn generated for recursive functions as well, and used in main fv for bindings.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1453
diff changeset
   169
  apply(simp_all add: eqvts)
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   170
  apply(simp add: alpha_gen)
1405
3e128904baba More tries about the proofs in trm5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1402
diff changeset
   171
  apply(clarify)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   172
  apply blast
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   173
done
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   174
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   175
lemma bv_list_rsp:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   176
  shows "x \<approx>l y \<Longrightarrow> rbv5 x = rbv5 y"
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   177
  apply(induct rule: alpha_rtrm5_alpha_rlts_alpha_rbv5.inducts(2))
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   178
  apply(simp_all)
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   179
  apply(clarify)
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   180
  apply simp
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   181
  done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   182
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   183
local_setup {* snd o Local_Theory.note ((@{binding alpha_dis}, []), (flat (map (distinct_rel @{context} @{thms alpha_rtrm5.cases alpha_rlts.cases alpha_rbv5.cases}) [(@{thms rtrm5.distinct}, @{term alpha_rtrm5}), (@{thms rlts.distinct}, @{term alpha_rlts}), (@{thms rlts.distinct}, @{term alpha_rbv5})]))) *}
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   184
print_theorems
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   185
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   186
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   187
lemma alpha_rbv_rsp_pre:
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   188
  "x \<approx>l y \<Longrightarrow> \<forall>z. alpha_rbv5 x z = alpha_rbv5 y z"
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   189
  apply (erule alpha_rtrm5_alpha_rlts_alpha_rbv5.inducts(2))
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   190
  apply (simp_all add: alpha_dis alpha5_inj)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   191
  apply clarify
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   192
  apply (case_tac [!] z)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   193
  apply (simp_all add: alpha_dis alpha5_inj)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   194
  apply clarify
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   195
  apply auto
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   196
  apply (meson alpha5_symp alpha5_transp)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   197
  apply (meson alpha5_symp alpha5_transp)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   198
  done
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   199
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   200
lemma alpha_rbv_rsp_pre2:
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   201
  "x \<approx>l y \<Longrightarrow> \<forall>z. alpha_rbv5 z x = alpha_rbv5 z y"
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   202
  apply (erule alpha_rtrm5_alpha_rlts_alpha_rbv5.inducts(2))
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   203
  apply (simp_all add: alpha_dis alpha5_inj)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   204
  apply clarify
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   205
  apply (case_tac [!] z)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   206
  apply (simp_all add: alpha_dis alpha5_inj)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   207
  apply clarify
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   208
  apply auto
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   209
  apply (meson alpha5_symp alpha5_transp)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   210
  apply (meson alpha5_symp alpha5_transp)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   211
  done
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   212
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   213
lemma [quot_respect]:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   214
  "(alpha_rlts ===> op =) fv_rlts fv_rlts"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   215
  "(alpha_rtrm5 ===> op =) fv_rtrm5 fv_rtrm5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   216
  "(alpha_rlts ===> op =) rbv5 rbv5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   217
  "(op = ===> alpha_rtrm5) rVr5 rVr5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   218
  "(alpha_rtrm5 ===> alpha_rtrm5 ===> alpha_rtrm5) rAp5 rAp5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   219
  "(alpha_rlts ===> alpha_rtrm5 ===> alpha_rtrm5) rLt5 rLt5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   220
  "(op = ===> alpha_rtrm5 ===> alpha_rlts ===> alpha_rlts) rLcons rLcons"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   221
  "(op = ===> alpha_rtrm5 ===> alpha_rtrm5) permute permute"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   222
  "(op = ===> alpha_rlts ===> alpha_rlts) permute permute"
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   223
  "(alpha_rlts ===> alpha_rlts ===> op =) alpha_rbv5 alpha_rbv5"
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   224
  apply (simp_all add: alpha5_inj alpha5_rfv alpha5_eqvt bv_list_rsp)
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   225
  apply (clarify)
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   226
  apply (rule_tac x="0" in exI)
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   227
  apply (simp add: fresh_star_def fresh_zero_perm alpha_gen alpha5_rfv)
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   228
  apply clarify
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   229
  apply (simp add: alpha_rbv_rsp_pre2)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   230
  apply (simp add: alpha_rbv_rsp_pre)
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   231
done
1405
3e128904baba More tries about the proofs in trm5
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1402
diff changeset
   232
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   233
lemma
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   234
  shows "(alpha_rlts ===> op =) rbv5 rbv5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   235
  by (simp add: bv_list_rsp)
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   236
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   237
lemmas trm5_lts_inducts = rtrm5_rlts.inducts[quot_lifted]
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   238
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   239
instantiation trm5 and lts :: pt
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   240
begin
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   241
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   242
quotient_definition
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   243
  "permute_trm5 :: perm \<Rightarrow> trm5 \<Rightarrow> trm5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   244
is
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   245
  "permute :: perm \<Rightarrow> rtrm5 \<Rightarrow> rtrm5"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   246
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   247
quotient_definition
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   248
  "permute_lts :: perm \<Rightarrow> lts \<Rightarrow> lts"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   249
is
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   250
  "permute :: perm \<Rightarrow> rlts \<Rightarrow> rlts"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   251
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   252
instance by default
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   253
  (simp_all add: permute_rtrm5_permute_rlts_zero[quot_lifted] permute_rtrm5_permute_rlts_append[quot_lifted])
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   254
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   255
end
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   256
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   257
lemmas permute_trm5_lts = permute_rtrm5_permute_rlts.simps[quot_lifted]
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   258
lemmas bv5[simp] = rbv5.simps[quot_lifted]
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   259
lemmas fv_trm5_lts[simp] = fv_rtrm5_fv_rlts.simps[quot_lifted]
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   260
lemmas alpha5_INJ = alpha5_inj[unfolded alpha_gen2, unfolded alpha_gen, quot_lifted, folded alpha_gen2, folded alpha_gen]
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   261
lemmas alpha5_DIS = alpha_dis[quot_lifted]
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   262
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   263
(* why is this not in Isabelle? *)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   264
lemma set_sub: "{a, b} - {b} = {a} - {b}"
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   265
by auto
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   266
1458
9cb619aa933c Alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1456
diff changeset
   267
lemma lets_bla:
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   268
  "x \<noteq> z \<Longrightarrow> y \<noteq> z \<Longrightarrow> x \<noteq> y \<Longrightarrow>(Lt5 (Lcons x (Vr5 y) Lnil) (Vr5 x)) \<noteq> (Lt5 (Lcons x (Vr5 z) Lnil) (Vr5 x))"
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   269
apply (simp only: alpha5_INJ bv5)
1458
9cb619aa933c Alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1456
diff changeset
   270
apply simp
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   271
apply (rule allI)
1458
9cb619aa933c Alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1456
diff changeset
   272
apply (simp_all add: alpha_gen)
9cb619aa933c Alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1456
diff changeset
   273
apply (simp add: permute_trm5_lts fresh_star_def alpha5_INJ eqvts)
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   274
apply (rule impI)
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   275
apply (rule impI)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   276
apply (rule impI)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   277
apply (simp add: set_sub)
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   278
done
1458
9cb619aa933c Alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1456
diff changeset
   279
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   280
lemma lets_ok:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   281
  "(Lt5 (Lcons x (Vr5 x) Lnil) (Vr5 x)) = (Lt5 (Lcons y (Vr5 y) Lnil) (Vr5 y))"
1454
7c8cd6eae8e2 FV_bn generated for recursive functions as well, and used in main fv for bindings.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1453
diff changeset
   282
thm alpha5_INJ
7c8cd6eae8e2 FV_bn generated for recursive functions as well, and used in main fv for bindings.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1453
diff changeset
   283
apply (simp only: alpha5_INJ)
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   284
apply (rule_tac x="(x \<leftrightarrow> y)" in exI)
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   285
apply (simp_all add: alpha_gen)
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   286
apply (simp add: permute_trm5_lts fresh_star_def)
1474
8a03753e0e02 Finished all proofs in Term5 and Term5n.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1464
diff changeset
   287
apply (simp add: eqvts)
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   288
done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   289
1286
87894b5156f4 Example that shows that current alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1277
diff changeset
   290
lemma lets_ok3:
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   291
  "x \<noteq> y \<Longrightarrow>
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   292
   (Lt5 (Lcons x (Ap5 (Vr5 y) (Vr5 x)) (Lcons y (Vr5 y) Lnil)) (Ap5 (Vr5 x) (Vr5 y))) \<noteq>
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   293
   (Lt5 (Lcons y (Ap5 (Vr5 x) (Vr5 y)) (Lcons x (Vr5 x) Lnil)) (Ap5 (Vr5 x) (Vr5 y)))"
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   294
apply (simp add: permute_trm5_lts alpha_gen alpha5_INJ)
1286
87894b5156f4 Example that shows that current alpha is wrong.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1277
diff changeset
   295
done
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   296
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   297
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   298
lemma lets_not_ok1:
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   299
  "x \<noteq> y \<Longrightarrow>
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   300
   (Lt5 (Lcons x (Vr5 x) (Lcons y (Vr5 y) Lnil)) (Ap5 (Vr5 x) (Vr5 y))) \<noteq>
1391
ebfbcadeac5e Testing equalities in trm5, all seems good.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1288
diff changeset
   301
   (Lt5 (Lcons y (Vr5 x) (Lcons x (Vr5 y) Lnil)) (Ap5 (Vr5 x) (Vr5 y)))"
1288
0203cd5cfd6c The new alpha-equivalence and testing in Trm2 and Trm5.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1287
diff changeset
   302
apply (simp add: alpha5_INJ alpha_gen)
1462
7c59dd8e5435 The old recursive alpha works fine.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1458
diff changeset
   303
apply (simp add: permute_trm5_lts eqvts)
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   304
apply (simp add: alpha5_INJ)
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   305
done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   306
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   307
lemma lets_nok:
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   308
  "x \<noteq> y \<Longrightarrow> x \<noteq> z \<Longrightarrow> z \<noteq> y \<Longrightarrow>
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   309
   (Lt5 (Lcons x (Ap5 (Vr5 z) (Vr5 z)) (Lcons y (Vr5 z) Lnil)) (Ap5 (Vr5 x) (Vr5 y))) \<noteq>
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   310
   (Lt5 (Lcons y (Vr5 z) (Lcons x (Ap5 (Vr5 z) (Vr5 z)) Lnil)) (Ap5 (Vr5 x) (Vr5 y)))"
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   311
apply (simp only: alpha5_INJ(3) alpha5_INJ(5) alpha_gen permute_trm5_lts fresh_star_def)
1464
1850361efb8f Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 1462
diff changeset
   312
apply (simp add: alpha5_DIS alpha5_INJ permute_trm5_lts)
1270
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   313
done
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   314
8c3cf9f4f5f2 Split Terms into separate files and add them to tests.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff changeset
   315
end