src/HOL/Nominal/Examples/SN.thy
changeset 29097 68245155eb58
parent 27272 75b251e9cdb7
child 32960 69916a850301
--- a/src/HOL/Nominal/Examples/SN.thy	Fri Dec 12 12:14:02 2008 +0100
+++ b/src/HOL/Nominal/Examples/SN.thy	Sat Dec 13 13:24:45 2008 +0100
@@ -1,5 +1,3 @@
-(* $Id$ *)
-
 theory SN
   imports Lam_Funs
 begin
@@ -228,12 +226,11 @@
 
 section {* Candidates *}
 
-consts
+nominal_primrec
   RED :: "ty \<Rightarrow> lam set"
-
-nominal_primrec
+where
   "RED (TVar X) = {t. SN(t)}"
-  "RED (\<tau>\<rightarrow>\<sigma>) =   {t. \<forall>u. (u\<in>RED \<tau> \<longrightarrow> (App t u)\<in>RED \<sigma>)}"
+| "RED (\<tau>\<rightarrow>\<sigma>) =   {t. \<forall>u. (u\<in>RED \<tau> \<longrightarrow> (App t u)\<in>RED \<sigma>)}"
 by (rule TrueI)+
 
 text {* neutral terms *}
@@ -248,13 +245,12 @@
 where
   fst[intro!]:  "(App t s) \<guillemotright> t"
 
-consts
+nominal_primrec
   fst_app_aux::"lam\<Rightarrow>lam option"
-
-nominal_primrec
+where
   "fst_app_aux (Var a)     = None"
-  "fst_app_aux (App t1 t2) = Some t1"
-  "fst_app_aux (Lam [x].t) = None"
+| "fst_app_aux (App t1 t2) = Some t1"
+| "fst_app_aux (Lam [x].t) = None"
 apply(finite_guess)+
 apply(rule TrueI)+
 apply(simp add: fresh_none)