src/HOL/Bali/State.thy
changeset 61424 c3658c18b7bc
parent 59807 22bc39064290
child 62042 6c6ccf573479
--- a/src/HOL/Bali/State.thy	Tue Oct 13 09:21:14 2015 +0200
+++ b/src/HOL/Bali/State.thy	Tue Oct 13 09:21:15 2015 +0200
@@ -143,7 +143,7 @@
 definition
   fields_table :: "prog \<Rightarrow> qtname \<Rightarrow> (fspec \<Rightarrow> field \<Rightarrow> bool)  \<Rightarrow> (fspec, ty) table" where
   "fields_table G C P =
-    map_option type \<circ> table_of (filter (split P) (DeclConcepts.fields G C))"
+    map_option type \<circ> table_of (filter (case_prod P) (DeclConcepts.fields G C))"
 
 lemma fields_table_SomeI: 
 "\<lbrakk>table_of (DeclConcepts.fields G C) n = Some f; P n f\<rbrakk>