diff -r 59b937edcff8 -r 4ec8e654112f src/HOL/Codegenerator_Test/Code_Lazy_Test.thy --- a/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Thu Jun 26 17:30:33 2025 +0200 +++ b/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Thu Jun 26 17:25:29 2025 +0200 @@ -112,7 +112,6 @@ definition f1 :: "bool \ bool \ bool \ nat llist \ unit" where "f1 _ _ _ _ = ()" -declare [[code drop: f1]] lemma f1_code1 [code]: "f1 b c d ns = Code.abort (STR ''4'') (\_. ())" "f1 b c True \<^bold>[n, m\<^bold>] = Code.abort (STR ''3'') (\_. ())" @@ -167,7 +166,6 @@ definition f2 :: "nat llist llist list \ unit" where "f2 _ = ()" -declare [[code drop: f2]] lemma f2_code1 [code]: "f2 xs = Code.abort (STR ''a'') (\_. ())" "f2 [\<^bold>[\<^bold>[\<^bold>]\<^bold>]] = ()" @@ -182,7 +180,6 @@ definition f3 :: "nat set llist \ unit" where "f3 _ = ()" -declare [[code drop: f3]] lemma f3_code1 [code]: "f3 \<^bold>[\<^bold>] = ()" "f3 \<^bold>[A\<^bold>] = ()"